src/ZF/Constructible/L_axioms.thy
changeset 29223 e09c53289830
parent 21404 eb85850d3eb7
child 30729 461ee3e49ad3
--- a/src/ZF/Constructible/L_axioms.thy	Wed Dec 10 17:19:25 2008 +0100
+++ b/src/ZF/Constructible/L_axioms.thy	Thu Dec 11 18:30:26 2008 +0100
@@ -1,5 +1,4 @@
 (*  Title:      ZF/Constructible/L_axioms.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
 *)
 
@@ -100,7 +99,7 @@
   apply (rule L_nat)
   done
 
-interpretation M_trivial ["L"] by (rule M_trivial_L)
+interpretation L: M_trivial L by (rule M_trivial_L)
 
 (* Replaces the following declarations...
 lemmas rall_abs = M_trivial.rall_abs [OF M_trivial_L]