Skip to content

Commit

Permalink
Fix a Moscow ML compilation error from recent changes
Browse files Browse the repository at this point in the history
  • Loading branch information
mn200 committed Jan 23, 2025
1 parent 8f3db54 commit 6c4ef89
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/portableML/rawtheory/RawTheoryReader.sml
Original file line number Diff line number Diff line change
Expand Up @@ -94,9 +94,9 @@ fun raw_term_decode s =
decoding raw theorems
---------------------------------------------------------------------- *)

fun decclass 0 = DB_dtype.Axm
| decclass 1 = DB_dtype.Def
| decclass 2 = DB_dtype.Thm
fun decclass 0 = Axm
| decclass 1 = Def
| decclass 2 = Thm
| decclass i = raise TheoryReader ("Bad theorem class: "^Int.toString i)

val dep_decode : int raw_dep decoder = let
Expand Down

0 comments on commit 6c4ef89

Please sign in to comment.