src/Pure/Isar/proof_context.ML
changeset 47247 23654b331d5c
parent 47005 421760a1efe7
child 47275 fc95b8b6c260
--- a/src/Pure/Isar/proof_context.ML	Sun Apr 01 15:23:43 2012 +0200
+++ b/src/Pure/Isar/proof_context.ML	Sun Apr 01 18:01:19 2012 +0200
@@ -136,9 +136,9 @@
   val get_case: Proof.context -> string -> binding option list -> Rule_Cases.T
   val type_notation: bool -> Syntax.mode -> (typ * mixfix) list -> Proof.context -> Proof.context
   val notation: bool -> Syntax.mode -> (term * mixfix) list -> Proof.context -> Proof.context
-  val target_type_notation: bool -> Syntax.mode -> (typ * mixfix) list -> morphism ->
+  val generic_type_notation: bool -> Syntax.mode -> (typ * mixfix) list -> morphism ->
     Context.generic -> Context.generic
-  val target_notation: bool -> Syntax.mode -> (term * mixfix) list -> morphism ->
+  val generic_notation: bool -> Syntax.mode -> (term * mixfix) list -> morphism ->
     Context.generic -> Context.generic
   val class_alias: binding -> class -> Proof.context -> Proof.context
   val type_alias: binding -> string -> Proof.context -> Proof.context
@@ -970,7 +970,7 @@
 val type_notation = gen_notation (K type_syntax);
 val notation = gen_notation const_syntax;
 
-fun target_type_notation add mode args phi =
+fun generic_type_notation add mode args phi =
   let
     val args' = args |> map_filter (fn (T, mx) =>
       let
@@ -979,7 +979,7 @@
       in if similar then SOME (T', mx) else NONE end);
   in Context.mapping (Sign.type_notation add mode args') (type_notation add mode args') end;
 
-fun target_notation add mode args phi =
+fun generic_notation add mode args phi =
   let
     val args' = args |> map_filter (fn (t, mx) =>
       let val t' = Morphism.term phi t