Import of AFP for Isabelle 2021.

This commit is contained in:
Achim D. Brucker 2021-02-27 16:34:10 +00:00
부모 2863b3552a
커밋 1f29340b1b
5개의 변경된 파일7개의 추가작업 그리고 12개의 파일을 삭제

파일 보기

@ -68,12 +68,10 @@ lemma mutex_not_gval:
apply simp
apply simp
apply simp
apply (case_tac "s v")
apply (case_tac "s v'")
apply simp
apply (case_tac "s v'")
apply simp
apply simp
apply simp
apply (case_tac "s v")
apply (case_tac "s v")
apply (case_tac "s v'")
by auto

파일 보기

파일 보기

@ -1,5 +1,5 @@
\documentclass[10pt,DIV16,a4paper,abstract=true,twoside=semi,openright]{scrreprt}
\usepackage[USenglish]{babel}
\usepackage[english]{babel}
\usepackage[numbers, sort&compress]{natbib}
\usepackage{isabelle,isabellesym}
\usepackage{booktabs}
@ -22,8 +22,6 @@
\begingroup%
\def\isacharunderscore{\textunderscore}%
\section{#1 (\thy)}%
\def\isacharunderscore{-}%
\expandafter\label{sec:\isabellecontext}%
\endgroup%
}

파일 보기

@ -1,5 +1,5 @@
subsection{*Example*}
text{*This theory shows how contexts can be used to prove transition subsumption.*}
subsection\<open>Example\<close>
text\<open>This theory shows how contexts can be used to prove transition subsumption.\<close>
theory Drinks_Subsumption
imports "Extended_Finite_State_Machine_Inference.Subsumption" "Extended_Finite_State_Machines.Drinks_Machine_2"
begin
@ -74,7 +74,6 @@ next
apply clarify
apply (simp add: in_possible_steps[symmetric])
apply (simp add: drinks2_def)
apply clarsimp
apply (simp add: drinks2_def[symmetric])
apply (simp add: select_def can_take apply_updates_def)
using no_change_1_1 by fastforce

파일 보기

@ -704,7 +704,7 @@ next
apply (induct a)
apply simp
apply simp
subgoal for _ x2 i ia
subgoal for x2 i ia
apply (case_tac x2)
apply (rule_tac x="list_update i ia x1" in exI)
apply (simp add: apply_guards_cons unconstrained_input filter_empty_conv)