Skip to content

Commit

Permalink
Modernise a theorem's syntax
Browse files Browse the repository at this point in the history
  • Loading branch information
mn200 committed Feb 3, 2023
1 parent fbf6a07 commit ff6e145
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/coalgebras/llistScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -744,10 +744,10 @@ val _ = computeLib.add_persistent_funs ["LAPPEND"]

(* properties of map and append *)

val LMAP_APPEND = store_thm(
"LMAP_APPEND",
``!f ll1 ll2. LMAP f (LAPPEND ll1 ll2) =
LAPPEND (LMAP f ll1) (LMAP f ll2)``,
Theorem LMAP_APPEND:
!f ll1 ll2.
LMAP f (LAPPEND ll1 ll2) = LAPPEND (LMAP f ll1) (LMAP f ll2)
Proof
REPEAT GEN_TAC THEN ONCE_REWRITE_TAC [LLIST_BISIMULATION0] THEN
Q.EXISTS_TAC `\ll1 ll2. ?x y. (ll1 = LMAP f (LAPPEND x y)) /\
(ll2 = LAPPEND (LMAP f x) (LMAP f y))` THEN
Expand Down

0 comments on commit ff6e145

Please sign in to comment.