src/HOL/Statespace/state_space.ML
changeset 74588 3cc363e8bfb2
parent 74586 5ac762b53119
child 78028 0ee49c509fea
equal deleted inserted replaced
74587:ebb0b15c66e1 74588:3cc363e8bfb2
     1 (*  Title:      HOL/Statespace/state_space.ML
     1 (*  Title:      HOL/Statespace/state_space.ML
     2     Author:     Norbert Schirmer, TU Muenchen
     2     Author:     Norbert Schirmer, TU Muenchen, 2007
       
     3     Author:     Norbert Schirmer, Apple, 2021
     3 *)
     4 *)
     4 
     5 
     5 signature STATE_SPACE =
     6 signature STATE_SPACE =
     6 sig
     7 sig
     7   val distinct_compsN : string
     8   val distinct_compsN : string
   657         Syntax.free (project_name T) $ Syntax.free n $ s
   658         Syntax.free (project_name T) $ Syntax.free n $ s
   658   | NONE =>
   659   | NONE =>
   659       if get_silent (Context.Proof ctxt)
   660       if get_silent (Context.Proof ctxt)
   660       then Syntax.const \<^const_name>\<open>StateFun.lookup\<close> $
   661       then Syntax.const \<^const_name>\<open>StateFun.lookup\<close> $
   661         Syntax.const \<^const_syntax>\<open>undefined\<close> $ Syntax.free n $ s
   662         Syntax.const \<^const_syntax>\<open>undefined\<close> $ Syntax.free n $ s
   662       else (trace_name_space_data (Context.Proof ctxt);
   663       else raise TERM ("StateSpace.gen_lookup_tr: component " ^ quote n ^ " not defined", []));
   663             raise TERM ("StateSpace.gen_lookup_tr: component " ^ quote n ^ " not defined", [])));
       
   664 
   664 
   665 fun lookup_tr ctxt [s, x] =
   665 fun lookup_tr ctxt [s, x] =
   666   (case Term_Position.strip_positions x of
   666   (case Term_Position.strip_positions x of
   667     Free (n,_) => gen_lookup_tr ctxt s n
   667     Free (n,_) => gen_lookup_tr ctxt s n
   668   | _ => raise Match);
   668   | _ => raise Match);