fixed type alias in signature;
authorwenzelm
Fri, 07 Sep 2007 20:40:08 +0200
changeset 24554 e9edafca311c
parent 24553 9b19da7b2b08
child 24555 ea220faa69e7
fixed type alias in signature;
src/Pure/Isar/local_theory.ML
--- a/src/Pure/Isar/local_theory.ML	Fri Sep 07 17:56:03 2007 +0200
+++ b/src/Pure/Isar/local_theory.ML	Fri Sep 07 20:40:08 2007 +0200
@@ -37,7 +37,7 @@
   val def: string -> (bstring * mixfix) * ((bstring * Attrib.src list) * term) ->
     local_theory -> (term * (bstring * thm)) * local_theory
   val note: string -> (bstring * Attrib.src list) * thm list ->
-    local_theory -> (bstring * thm list) * Proof.context
+    local_theory -> (bstring * thm list) * local_theory
   val notation: Syntax.mode -> (term * mixfix) list -> local_theory -> local_theory
   val target_morphism: local_theory -> morphism
   val target_naming: local_theory -> NameSpace.naming